// This prints the left floatting menu
Dedukti    Load Matita      Load Coq         Load Lean        Load PVS         Load OpenTheory Load
Dedukti-jumb

Theorem

fermat.prime_to_not_divides_fact

Statement

∀ p, prime p ⇒ ∀ n, n < p ⇒ ¬(p | (!n))

Main Dependencies
Theory

Coq-Jumb
Statement

Theorem prime_to_not_divides_fact : forall (p:nat.nat), (primes.prime p) -> forall (n:nat.nat), (nat.lt n p) -> connectives.Not (primes.divides p (fact.fact n)).



Matita-Jumb
Statement

theorem prime_to_not_divides_fact : \forall (p:nat). ((prime) p) -> \forall (n:nat). ((lt) n p) -> (Not) ((divides) p ((fact) n)).



Lean-jumb
Statement

theorem prime_to_not_divides_fact : forall (p:nat.nat) , (((primes.prime) ) (p)) -> forall (n:nat.nat) , ((((nat.lt_) ) (n)) (p)) -> ((connectives.Not) ) ((((primes.divides) ) (p)) (((fact.fact) ) (n))).



PVS-jumb

Statement

prime_to_not_divides_fact : LEMMA (FORALL(p:nat_sttfa_th.sttfa_nat):(primes_sttfa_th.prime(p) => (FORALL(n:nat_sttfa_th.sttfa_nat):(nat_sttfa_th.lt(n)(p) => connectives_sttfa_th.sttfa_Not(primes_sttfa_th.sttfa_divides(p)(fact_sttfa_th.sttfa_fact(n)))))))



OpenTheory

Printing for OpenTheory is not working at the moment.