src/HOL/List.thy
changeset 62100 7a5754afe170
parent 62090 db9996a84166
parent 62093 bd73a2279fcd
child 62175 8ffc4d0e652d
equal deleted inserted replaced
62090:db9996a84166 62100:7a5754afe170
  5650 
  5650 
  5651 context ord
  5651 context ord
  5652 begin
  5652 begin
  5653 
  5653 
  5654 context
  5654 context
  5655   notes [[inductive_defs]]
  5655   notes [[inductive_internals]]
  5656 begin
  5656 begin
  5657 
  5657 
  5658 inductive lexordp :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool"
  5658 inductive lexordp :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool"
  5659 where
  5659 where
  5660   Nil: "lexordp [] (y # ys)"
  5660   Nil: "lexordp [] (y # ys)"