From 9058fb97426307536f56c3e7447be2f70798e081 Mon Sep 17 00:00:00 2001 From: herbelin Date: Sat, 29 Nov 2003 16:15:58 +0000 Subject: Deplacement des fichiers ancienne syntaxe dans theories7, contrib7 et states7 git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5026 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories7/Sets/Relations_3.v | 63 ++++++++++++++++++++++++++++++++++++++++++++ 1 file changed, 63 insertions(+) create mode 100755 theories7/Sets/Relations_3.v (limited to 'theories7/Sets/Relations_3.v') diff --git a/theories7/Sets/Relations_3.v b/theories7/Sets/Relations_3.v new file mode 100755 index 000000000..90c055775 --- /dev/null +++ b/theories7/Sets/Relations_3.v @@ -0,0 +1,63 @@ +(***********************************************************************) +(* v * The Coq Proof Assistant / The Coq Development Team *) +(* U -> Prop := + [x,y: U] (EXT z | (Rstar U R x z) /\ (Rstar U R y z)). + + Definition locally_confluent : U -> Prop := + [x: U] (y,z: U) (R x y) -> (R x z) -> (coherent y z). + + Definition Locally_confluent : Prop := (x: U) (locally_confluent x). + + Definition confluent : U -> Prop := + [x: U] (y,z: U) (Rstar U R x y) -> (Rstar U R x z) -> (coherent y z). + + Definition Confluent : Prop := (x: U) (confluent x). + + Inductive noetherian : U -> Prop := + definition_of_noetherian: + (x: U) ((y: U) (R x y) -> (noetherian y)) -> (noetherian x). + + Definition Noetherian : Prop := (x: U) (noetherian x). + +End Relations_3. +Hints Unfold coherent : sets v62. +Hints Unfold locally_confluent : sets v62. +Hints Unfold confluent : sets v62. +Hints Unfold Confluent : sets v62. +Hints Resolve definition_of_noetherian : sets v62. +Hints Unfold Noetherian : sets v62. + + -- cgit v1.2.3