src/HOL/Codegenerator_Test/Candidates.thy
changeset 41884 335895ffbd94
parent 37695 71e84a203c19
child 49077 154f25a162e3
equal deleted inserted replaced
41883:392364739e5d 41884:335895ffbd94
     5 
     5 
     6 theory Candidates
     6 theory Candidates
     7 imports
     7 imports
     8   Complex_Main
     8   Complex_Main
     9   Library
     9   Library
    10   List_Prefix
    10   "~~/src/HOL/Library/List_Prefix"
    11   "~~/src/HOL/Number_Theory/Primes"
    11   "~~/src/HOL/Number_Theory/Primes"
    12   "~~/src/HOL/ex/Records"
    12   "~~/src/HOL/ex/Records"
    13 begin
    13 begin
    14 
    14 
    15 inductive sublist :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool" where
    15 inductive sublist :: "'a list \<Rightarrow> 'a list \<Rightarrow> bool" where