src/HOL/Library/Dense_Linear_Order.thy
changeset 26199 04817a8802f2
parent 26161 34cb0b457dcc
child 27368 9f90ac19e32b
equal deleted inserted replaced
26198:865bca530d4c 26199:04817a8802f2
   262   using gt_ex[of t] by auto
   262   using gt_ex[of t] by auto
   263 
   263 
   264 lemmas dlo_simps = order_refl less_irrefl not_less not_le exists_neq 
   264 lemmas dlo_simps = order_refl less_irrefl not_less not_le exists_neq 
   265   le_less neq_iff linear less_not_permute
   265   le_less neq_iff linear less_not_permute
   266 
   266 
   267 lemma axiom: "dense_linear_order (op \<le>) (op <)" by fact
   267 lemma axiom: "dense_linear_order (op \<le>) (op <)" by (rule dense_linear_order_axioms)
   268 lemma atoms:
   268 lemma atoms:
   269   includes meta_term_syntax
   269   includes meta_term_syntax
   270   shows "TERM (less :: 'a \<Rightarrow> _)"
   270   shows "TERM (less :: 'a \<Rightarrow> _)"
   271     and "TERM (less_eq :: 'a \<Rightarrow> _)"
   271     and "TERM (less_eq :: 'a \<Rightarrow> _)"
   272     and "TERM (op = :: 'a \<Rightarrow> _)" .
   272     and "TERM (op = :: 'a \<Rightarrow> _)" .
   498 
   498 
   499 lemmas nmi_thms = nmi_conj nmi_disj nmi_eq nmi_neq nmi_lt nmi_le nmi_gt nmi_ge nmi_P
   499 lemmas nmi_thms = nmi_conj nmi_disj nmi_eq nmi_neq nmi_lt nmi_le nmi_gt nmi_ge nmi_P
   500 lemmas npi_thms = npi_conj npi_disj npi_eq npi_neq npi_lt npi_le npi_gt npi_ge npi_P
   500 lemmas npi_thms = npi_conj npi_disj npi_eq npi_neq npi_lt npi_le npi_gt npi_ge npi_P
   501 lemmas lin_dense_thms = lin_dense_conj lin_dense_disj lin_dense_eq lin_dense_neq lin_dense_lt lin_dense_le lin_dense_gt lin_dense_ge lin_dense_P
   501 lemmas lin_dense_thms = lin_dense_conj lin_dense_disj lin_dense_eq lin_dense_neq lin_dense_lt lin_dense_le lin_dense_gt lin_dense_ge lin_dense_P
   502 
   502 
   503 lemma ferrack_axiom: "constr_dense_linear_order less_eq less between" by fact
   503 lemma ferrack_axiom: "constr_dense_linear_order less_eq less between"
       
   504   by (rule constr_dense_linear_order_axioms)
   504 lemma atoms:
   505 lemma atoms:
   505   includes meta_term_syntax
   506   includes meta_term_syntax
   506   shows "TERM (less :: 'a \<Rightarrow> _)"
   507   shows "TERM (less :: 'a \<Rightarrow> _)"
   507     and "TERM (less_eq :: 'a \<Rightarrow> _)"
   508     and "TERM (less_eq :: 'a \<Rightarrow> _)"
   508     and "TERM (op = :: 'a \<Rightarrow> _)" .
   509     and "TERM (op = :: 'a \<Rightarrow> _)" .