From 6b649aba925b6f7462da07599fe67ebb12a3460e Mon Sep 17 00:00:00 2001 From: Samuel Mimram Date: Wed, 28 Jul 2004 21:54:47 +0000 Subject: Imported Upstream version 8.0pl1 --- 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 00000000..092fc534 --- /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