src/HOL/BNF_Wellorder_Constructions.thy
changeset 63561 fba08009ff3e
parent 63092 a949b2a5f51d
child 67091 1393c2340eec
--- a/src/HOL/BNF_Wellorder_Constructions.thy	Thu Jul 28 20:39:51 2016 +0200
+++ b/src/HOL/BNF_Wellorder_Constructions.thy	Fri Jul 29 09:49:23 2016 +0200
@@ -36,6 +36,10 @@
 lemma Refl_Restr: "Refl r \<Longrightarrow> Refl(Restr r A)"
 unfolding refl_on_def Field_def by auto
 
+lemma linear_order_on_Restr:
+  "linear_order_on A r \<Longrightarrow> linear_order_on (A \<inter> above r x) (Restr r (above r x))"
+by(simp add: order_on_defs refl_on_def trans_def antisym_def total_on_def)(safe; blast)
+
 lemma antisym_Restr:
 "antisym r \<Longrightarrow> antisym(Restr r A)"
 unfolding antisym_def Field_def by auto